coq

    20Hitze

    5Antwort

    Kennt jemand Beispiele für die folgenden? Proof Entwicklungen über regular expressions (evtl. mit backreferences erweitert) in Beweisassistenten (wie Coq). Programme in abhängigen Sprachen (z. B. Agda

    2Hitze

    2Antwort

    Ich versuche Coq, aber ich bin mir nicht ganz sicher, was ich mache. Ist: Theorem new_theorem : forall x, P:Prop /\ Q:Prop Entspricht: ∀x (P(x) and Q(x)) Edit: Ich denke, sie sind.

    5Hitze

    1Antwort

    Ich habe die definierten induktiven Typen: Inductive InL (A:Type) (y:A) : list A -> Prop := | InHead : forall xs:list A, InL y (cons y xs) | InTail : forall (x:A) (xs:list A), InL y xs -> In