doc-src/IsarImplementation/Thy/Isar.thy
changeset 40149 4c35be108990
parent 40126 916cb4a28ffd
child 40800 330eb65c9469
equal deleted inserted replaced
40148:8728165d366e 40149:4c35be108990
   359   \cite{isabelle-isar-ref} which includes some abstract examples.
   359   \cite{isabelle-isar-ref} which includes some abstract examples.
   360 
   360 
   361   \medskip The following toy examples illustrate how the goal facts
   361   \medskip The following toy examples illustrate how the goal facts
   362   and state are passed to proof methods.  The pre-defined proof method
   362   and state are passed to proof methods.  The pre-defined proof method
   363   called ``@{method tactic}'' wraps ML source of type @{ML_type
   363   called ``@{method tactic}'' wraps ML source of type @{ML_type
   364   tactic} (abstracted over @{verbatim facts}).  This allows immediate
   364   tactic} (abstracted over @{ML_text facts}).  This allows immediate
   365   experimentation without parsing of concrete syntax. *}
   365   experimentation without parsing of concrete syntax. *}
   366 
   366 
   367 example_proof
   367 example_proof
   368   assume a: A and b: B
   368   assume a: A and b: B
   369 
   369 
   396   not used in this example.
   396   not used in this example.
   397 
   397 
   398   The @{ML Attrib.thms} parser produces a list of theorems from the
   398   The @{ML Attrib.thms} parser produces a list of theorems from the
   399   usual Isar syntax involving attribute expressions etc.\ (syntax
   399   usual Isar syntax involving attribute expressions etc.\ (syntax
   400   category @{syntax thmrefs}) \cite{isabelle-isar-ref}.  The resulting
   400   category @{syntax thmrefs}) \cite{isabelle-isar-ref}.  The resulting
   401   @{verbatim thms} are added to @{ML HOL_basic_ss} which already
   401   @{ML_text thms} are added to @{ML HOL_basic_ss} which already
   402   contains the basic Simplifier setup for HOL.
   402   contains the basic Simplifier setup for HOL.
   403 
   403 
   404   The tactic @{ML asm_full_simp_tac} is the one that is also used in
   404   The tactic @{ML asm_full_simp_tac} is the one that is also used in
   405   method @{method simp} by default.  The extra wrapping by the @{ML
   405   method @{method simp} by default.  The extra wrapping by the @{ML
   406   CHANGED} tactical ensures progress of simplification: identical goal
   406   CHANGED} tactical ensures progress of simplification: identical goal