doc-src/IsarRef/Thy/Generic.thy
changeset 47497 c78c6e1ec75d
parent 46706 877d57975427
child 47967 c422128d3889
equal deleted inserted replaced
47496:a43f207f216f 47497:c78c6e1ec75d
   127     @{attribute_def tagged} & : & @{text attribute} \\
   127     @{attribute_def tagged} & : & @{text attribute} \\
   128     @{attribute_def untagged} & : & @{text attribute} \\[0.5ex]
   128     @{attribute_def untagged} & : & @{text attribute} \\[0.5ex]
   129     @{attribute_def THEN} & : & @{text attribute} \\
   129     @{attribute_def THEN} & : & @{text attribute} \\
   130     @{attribute_def COMP} & : & @{text attribute} \\[0.5ex]
   130     @{attribute_def COMP} & : & @{text attribute} \\[0.5ex]
   131     @{attribute_def unfolded} & : & @{text attribute} \\
   131     @{attribute_def unfolded} & : & @{text attribute} \\
   132     @{attribute_def folded} & : & @{text attribute} \\[0.5ex]
   132     @{attribute_def folded} & : & @{text attribute} \\
       
   133     @{attribute_def abs_def} & : & @{text attribute} \\[0.5ex]
   133     @{attribute_def rotated} & : & @{text attribute} \\
   134     @{attribute_def rotated} & : & @{text attribute} \\
   134     @{attribute_def (Pure) elim_format} & : & @{text attribute} \\
   135     @{attribute_def (Pure) elim_format} & : & @{text attribute} \\
   135     @{attribute_def standard}@{text "\<^sup>*"} & : & @{text attribute} \\
   136     @{attribute_def standard}@{text "\<^sup>*"} & : & @{text attribute} \\
   136     @{attribute_def no_vars}@{text "\<^sup>*"} & : & @{text attribute} \\
   137     @{attribute_def no_vars}@{text "\<^sup>*"} & : & @{text attribute} \\
   137   \end{matharray}
   138   \end{matharray}
   164   @{ML_op "COMP"} in \cite{isabelle-implementation}).
   165   @{ML_op "COMP"} in \cite{isabelle-implementation}).
   165   
   166   
   166   \item @{attribute unfolded}~@{text "a\<^sub>1 \<dots> a\<^sub>n"} and @{attribute
   167   \item @{attribute unfolded}~@{text "a\<^sub>1 \<dots> a\<^sub>n"} and @{attribute
   167   folded}~@{text "a\<^sub>1 \<dots> a\<^sub>n"} expand and fold back again the given
   168   folded}~@{text "a\<^sub>1 \<dots> a\<^sub>n"} expand and fold back again the given
   168   definitions throughout a rule.
   169   definitions throughout a rule.
       
   170 
       
   171   \item @{attribute abs_def} turns an equation of the form @{prop "f x
       
   172   y \<equiv> t"} into @{prop "f \<equiv> \<lambda>x y. t"}, which ensures that @{method
       
   173   simp} or @{method unfold} steps always expand it.  This also works
       
   174   for object-logic equality.
   169 
   175 
   170   \item @{attribute rotated}~@{text n} rotate the premises of a
   176   \item @{attribute rotated}~@{text n} rotate the premises of a
   171   theorem by @{text n} (default 1).
   177   theorem by @{text n} (default 1).
   172 
   178 
   173   \item @{attribute (Pure) elim_format} turns a destruction rule into
   179   \item @{attribute (Pure) elim_format} turns a destruction rule into