# Script simulating a dialog between coqide and coqtop -ideslave
# Run it via fake_ide
#
# Bug 2082
# Broken due to proof engine rewriting
#
ADD { Variable A : Prop. }
ADD { Variable B : Prop. }
ADD { Axiom OR : A \/ B. }
ADD { Lemma MyLemma2 : True. }
ADD { proof. }
ADD { per cases of (A \/ B) by OR. }
ADD { suppose A. }
ADD { then (1 = 1). }
ADD there { then H1 : thesis. }
ADD here { thus thesis by H1. }
ADD { suppose B. }
QUERY { Show. }
EDIT_AT here
#
ADD { suppose B. }
#
EDIT_AT there
#
ADD { thus thesis by H1. }
ADD { suppose B. }
#
QUERY { Show. }
ADD { then (1 = 1). }
ADD { then H2 : thesis. }
ADD { thus thesis by H2. }
ADD { end cases. }
ADD { end proof. }
ADD { Qed. }