doc-src/ZF/FOL_examples.thy
changeset 16417 9bc16273c2d4
parent 14152 12f6f18e7afc
child 48517 0f8c8ac6cc0e
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     1 header{*Examples of Classical Reasoning*}
     1 header{*Examples of Classical Reasoning*}
     2 
     2 
     3 theory FOL_examples = FOL:
     3 theory FOL_examples imports FOL begin
     4 
     4 
     5 lemma "EX y. ALL x. P(y)-->P(x)"
     5 lemma "EX y. ALL x. P(y)-->P(x)"
     6   --{* @{subgoals[display,indent=0,margin=65]} *}
     6   --{* @{subgoals[display,indent=0,margin=65]} *}
     7 apply (rule exCI)
     7 apply (rule exCI)
     8   --{* @{subgoals[display,indent=0,margin=65]} *}
     8   --{* @{subgoals[display,indent=0,margin=65]} *}