Skip to content

Commit

Permalink
clean up
Browse files Browse the repository at this point in the history
  • Loading branch information
tomaz1502 committed Oct 24, 2023
1 parent 690be60 commit 34385c4
Showing 1 changed file with 0 additions and 8 deletions.
8 changes: 0 additions & 8 deletions Smt/Tactic/Cvc5Proof.lean
Original file line number Diff line number Diff line change
Expand Up @@ -135,11 +135,6 @@ def cvc5Proof4: Cvc5Proof := {
lastName := `pf
}

example (P Q : Prop) : Q → ¬ P ∨ Q := by
intro lean_a0
have lean_a1: ¬ P ∨ Q := scope (fun hp => lean_a0)
exact lean_a1

def cvc5Proof5: Cvc5Proof := {
steps := [ .intro `lean_a0
, .scope `lean_a1 "P" "Q" `hp `inner_pf
Expand Down Expand Up @@ -176,6 +171,3 @@ example (P Q : Prop) : Not (P → ((P → Q) → Q)) → False := by
example (P Q : Prop) : Q → ¬ P ∨ Q := by
test 5

/- intro lean_a0 -/
/- have lean_a1: ¬ P ∨ Q := scope (fun hp => lean_a0) -/
/- exact lean_a1 -/

0 comments on commit 34385c4

Please sign in to comment.