changeset 80914 | d97fdabd9e2b |
parent 74888 | 1c50ddcf6a01 |
--- a/src/HOL/Library/Rewrite.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Library/Rewrite.thy Fri Sep 20 19:51:08 2024 +0200 @@ -10,7 +10,7 @@ imports Main begin -consts rewrite_HOLE :: "'a::{}" ("\<hole>") +consts rewrite_HOLE :: "'a::{}" (\<open>\<hole>\<close>) lemma eta_expand: fixes f :: "'a::{} \<Rightarrow> 'b::{}"